src/HOLCF/Lift1.ML
author oheimb
Wed, 18 Dec 1996 15:16:13 +0100
changeset 2445 51993fea433f
parent 2357 dd2e5e655fd2
child 2640 ee4dfce170a0
permissions -rw-r--r--
removed Holcfb.thy and Holcfb.ML, moving classical3 to HOL.ML as classical2

(*  Title:      HOLCF/Lift1.ML
    ID:         $Id$
    Author:     Olaf Mueller, Robert Sandner
    Copyright   1996 Technische Universitaet Muenchen

Theorems for Lift1.thy
*)


open Lift1;

(* ------------------------------------------------------------------------ *)
(* less_lift is a partial order on type 'a -> 'b                            *)
(* ------------------------------------------------------------------------ *)

goalw Lift1.thy [less_lift_def] "less_lift x x";
by (fast_tac HOL_cs 1);
qed"refl_less_lift";

goalw Lift1.thy [less_lift_def] 
  "less_lift x1 x2 & less_lift x2 x1 --> x1 = x2";
by (fast_tac HOL_cs 1);
qed"antisym_less_lift";

goalw Lift1.thy [less_lift_def] 
  "less_lift x1 x2 & less_lift x2 x3 --> less_lift x1 x3";
by (fast_tac HOL_cs 1);
qed"trans_less_lift";