src/HOLCF/FOCUS/FOCUS.ML
author kleing
Mon, 21 Jun 2004 10:25:57 +0200
changeset 14981 e73f8140af78
parent 12039 ef2a6fdd3564
child 15188 9d57263faf9e
permissions -rw-r--r--
Merged in license change from Isabelle2004

(*  Title: 	HOLCF/FOCUS/FOCUS.ML
    ID:         $Id$
    Author: 	David von Oheimb, TU Muenchen
*)

val ex_eqI = prove_goal thy "? xx. x = xx" (K [Auto_tac]);
val ex2_eqI = prove_goal thy "? xx yy. x = xx & y = yy" (K [Auto_tac]);
val eq_UU_symf = prove_goal thy "(UU = f x) = (f x = UU)" (K [Auto_tac]);

AddSIs [ex_eqI, ex2_eqI];
Addsimps[eq_UU_symf];
Goal "(#x ~= 0) = (? a y. x = a~> y)";
by (simp_tac (simpset() addsimps [slen_empty_eq, fstream_exhaust_eq]) 1);
qed "fstream_exhaust_slen_eq";

Addsimps[slen_less_1_eq, fstream_exhaust_slen_eq,
		   slen_fscons_eq, slen_fscons_less_eq];
Addsimps[thm "Suc_ile_eq"];
AddEs  [strictI];