Skip to content
Snippets Groups Projects
Commit 8bd02d0f authored by Ralf Jung's avatar Ralf Jung
Browse files

compile again

parent cf4310ed
No related branches found
No related tags found
No related merge requests found
(** This file provides the proof that CBUlt, the category of complete, (** This file provides the proof that CBUlt, the category of complete,
bisected, ultrametric spaces, forms an M-category. *) bisected, ultrametric spaces, forms an M-category. *)
Require Import MetricCore. Require Import CSetoid Constr.
Require Import MetricRec. Require Import MetricCore MetricRec.
Module CBUlt <: MCat. Module CBUlt <: MCat.
Local Open Scope cat_scope. Local Open Scope cat_scope.
......
...@@ -6,16 +6,9 @@ ...@@ -6,16 +6,9 @@
- an extension operation on the space Tᵏ, for k ∈ nat, as a - an extension operation on the space Tᵏ, for k ∈ nat, as a
non-expansive morphism. *) non-expansive morphism. *)
Require Export UPred. Require Import UPred.
Require Import MetricCore. Require Import MetricCore.
Require Import Arith. Require Fin.
Module NatDec.
Definition U := nat.
Definition eq_dec := eq_nat_dec.
End NatDec.
Module D := Coq.Logic.Eqdep_dec.DecidableEqDep(NatDec).
Section Halving. Section Halving.
Context (T : cmtyp). Context (T : cmtyp).
...@@ -174,8 +167,6 @@ Section EvaluationClosure. ...@@ -174,8 +167,6 @@ Section EvaluationClosure.
End EvaluationClosure. End EvaluationClosure.
Require Fin.
Definition transfer {A} {T : A -> Type} {x y : A} (EQ : x = y) (t : T x) : T y := Definition transfer {A} {T : A -> Type} {x y : A} (EQ : x = y) (t : T x) : T y :=
eq_rect x T t y EQ. eq_rect x T t y EQ.
......
...@@ -1001,3 +1001,11 @@ Section Option. ...@@ -1001,3 +1001,11 @@ Section Option.
End Option. End Option.
Arguments dist {_ _ _} _ _ _ /. Arguments dist {_ _ _} _ _ _ /.
(* We have several users of this, so deifne it centrally *)
Module NatDec.
Definition U := nat.
Definition eq_dec := eq_nat_dec.
End NatDec.
Module D := Coq.Logic.Eqdep_dec.DecidableEqDep(NatDec).
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment