aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--Makefile.common2
-rw-r--r--tactics/class_setoid.ml48
-rw-r--r--theories/Classes/SetoidClass.v (renamed from theories/Classes/Setoid.v)0
-rw-r--r--theories/Classes/SetoidTactics.v2
4 files changed, 6 insertions, 6 deletions
diff --git a/Makefile.common b/Makefile.common
index 84a15bf83..a8801f3df 100644
--- a/Makefile.common
+++ b/Makefile.common
@@ -706,7 +706,7 @@ SETOIDSVO:= theories/Setoids/Setoid_tac.vo theories/Setoids/Setoid_Prop.vo theor
UNICODEVO:= theories/Unicode/Utf8.vo
-CLASSESVO:= theories/Classes/Init.vo theories/Classes/Setoid.vo theories/Classes/SetoidTactics.v
+CLASSESVO:= theories/Classes/Init.vo theories/Classes/SetoidClass.vo theories/Classes/SetoidTactics.v
THEORIESVO:=\
$(INITVO) $(LOGICVO) $(ARITHVO) $(BOOLVO) $(NARITHVO) $(ZARITHVO) \
diff --git a/tactics/class_setoid.ml4 b/tactics/class_setoid.ml4
index 0c8bdd298..9111ba97e 100644
--- a/tactics/class_setoid.ml4
+++ b/tactics/class_setoid.ml4
@@ -57,10 +57,10 @@ let coq_proj1 = lazy(gen_constant ["Init"; "Logic"] "proj1")
let coq_proj2 = lazy(gen_constant ["Init"; "Logic"] "proj2")
let iff = lazy (gen_constant ["Init"; "Logic"] "iff")
-let iff_setoid = lazy (gen_constant ["Classes"; "Setoid"] "iff_setoid")
-let setoid_equiv = lazy (gen_constant ["Classes"; "Setoid"] "equiv")
-let setoid_morphism = lazy (gen_constant ["Classes"; "Setoid"] "setoid_morphism")
-let setoid_refl_proj = lazy (gen_constant ["Classes"; "Setoid"] "equiv_refl")
+let iff_setoid = lazy (gen_constant ["Classes"; "SetoidClass"] "iff_setoid")
+let setoid_equiv = lazy (gen_constant ["Classes"; "SetoidClass"] "equiv")
+let setoid_morphism = lazy (gen_constant ["Classes"; "SetoidClass"] "setoid_morphism")
+let setoid_refl_proj = lazy (gen_constant ["Classes"; "SetoidClass"] "equiv_refl")
let arrow_morphism a b =
mkLambda (Name (id_of_string "A"), a,
diff --git a/theories/Classes/Setoid.v b/theories/Classes/SetoidClass.v
index 915a7a944..915a7a944 100644
--- a/theories/Classes/Setoid.v
+++ b/theories/Classes/SetoidClass.v
diff --git a/theories/Classes/SetoidTactics.v b/theories/Classes/SetoidTactics.v
index 8e037db1a..4832f1d72 100644
--- a/theories/Classes/SetoidTactics.v
+++ b/theories/Classes/SetoidTactics.v
@@ -19,7 +19,7 @@ Require Import Coq.Program.Program.
Set Implicit Arguments.
Unset Strict Implicit.
-Require Export Coq.Classes.Setoid.
+Require Export Coq.Classes.SetoidClass.
Ltac rew H := clrewrite H.