# HG changeset patch # User wenzelm # Date 1444488043 -7200 # Node ID 6762c84451385086855dd38354d804258b665176 # Parent efac889fccbcfa34f01aa605a92635382fe1d87b use Isabelle symbols by default; diff -r efac889fccbc -r 6762c8445138 src/HOL/Library/Rewrite.thy --- a/src/HOL/Library/Rewrite.thy Sat Oct 10 16:26:23 2015 +0200 +++ b/src/HOL/Library/Rewrite.thy Sat Oct 10 16:40:43 2015 +0200 @@ -8,9 +8,7 @@ imports Main begin -consts rewrite_HOLE :: "'a::{}" -notation rewrite_HOLE ("HOLE") -notation rewrite_HOLE ("\") +consts rewrite_HOLE :: "'a::{}" ("\") lemma eta_expand: fixes f :: "'a::{} \ 'b::{}" @@ -25,7 +23,8 @@ done lemma imp_cong_eq: - "(PROP A \ (PROP B \ PROP C) \ (PROP B' \ PROP C')) \ ((PROP B \ PROP A \ PROP C) \ (PROP B' \ PROP A \ PROP C'))" + "(PROP A \ (PROP B \ PROP C) \ (PROP B' \ PROP C')) \ + ((PROP B \ PROP A \ PROP C) \ (PROP B' \ PROP A \ PROP C'))" apply (intro Pure.equal_intr_rule) apply (drule (1) cut_rl; drule Pure.equal_elim_rule1 Pure.equal_elim_rule2; assumption)+ apply (drule Pure.equal_elim_rule1 Pure.equal_elim_rule2; assumption)+