From 1eac679a065d9b161004fa4da881fdd734531693 Mon Sep 17 00:00:00 2001 From: notin Date: Thu, 16 Aug 2007 14:52:49 +0000 Subject: Correction du bug #1322 git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10077 85f007b7-540e-0410-9357-904b9bb8a0f7 --- test-suite/bugs/closed/1322.v | 24 ++++++++++++++++++++++++ 1 file changed, 24 insertions(+) create mode 100644 test-suite/bugs/closed/1322.v (limited to 'test-suite/bugs') diff --git a/test-suite/bugs/closed/1322.v b/test-suite/bugs/closed/1322.v new file mode 100644 index 000000000..01c06f2c4 --- /dev/null +++ b/test-suite/bugs/closed/1322.v @@ -0,0 +1,24 @@ +Require Import Setoid. + +Section transition_gen. + +Variable I : Type. +Variable I_eq :I -> I -> Prop. +Variable I_eq_equiv : Setoid_Theory I I_eq. + +(* Add Relation I I_eq + reflexivity proved by I_eq_equiv.(Seq_refl I I_eq) + symmetry proved by I_eq_equiv.(Seq_sym I I_eq) + transitivity proved by I_eq_equiv.(Seq_trans I I_eq) +as I_eq_relation. *) + +Add Setoid I I_eq I_eq_equiv as I_with_eq. + +Variable F : I -> Type. +Variable F_morphism : forall i j, I_eq i j -> F i = F j. + + +Add Morphism F with signature I_eq ==> eq as F_morphism2. +Admitted. + +End transition_gen. -- cgit v1.2.3