Lvc.Infra.Indexwise

Require Import Arith Coq.Lists.List Setoid Coq.Lists.SetoidList Omega Containers.OrderedTypeEx.
Require Export Infra.Option EqDec AutoIndTac Get.

Set Implicit Arguments.

Definition indexwise_R {A} {B} (R:ABProp) LA LB :=
n a b, get LA n aget LB n bR a b.

Definition indexwise_R_dec {A} {B} {R:ABProp} (Rdec:( a b, Computable (R a b))) LA LB
      : Computable (indexwise_R R LA LB) .
Defined.

Definition indexwise_R_dec´ {A} {B} {R:ABProp} LA LB (Rdec:( n a b, get LA n aget LB n bComputable (R a b)))
      : Computable (indexwise_R R LA LB).
Defined.